You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
import tactic
example (X : Type) (p : X → Prop) : (∃ x, p x) ↔ ¬ (∀ x, ¬ p x) :=
begin
library_search -- avoid smileys if you want to use "try this" :-)endexample (X : Type) (p : X → Prop) : (∃ x, p x) ↔ ¬ (∀ x, ¬ p x) :=
begin
library_search -- and frownies are even worse :-(end
Clicking on the "Try this:" code doesn't work, because the system gets confused by the brackets (in the first case the comment is deleted apart from the bracket; in the second case end gets deleted too). In practice I guess one isn't going to write anything after library_search usually -- the only reason I ran into this was because I was documenting something for a beginner.
Clicking on the "Try this:" code doesn't work, because the system gets confused by the brackets (in the first case the comment is deleted apart from the bracket; in the second case
end
gets deleted too). In practice I guess one isn't going to write anything after library_search usually -- the only reason I ran into this was because I was documenting something for a beginner.Originally opened by @kbuzzard as leanprover-community/mathlib3#5051
The text was updated successfully, but these errors were encountered: