c133d26505
Unresolved placeholders were not being reported
7 lines
185 B
Text
7 lines
185 B
Text
example (a b : Prop) : a ∧ b → b ∧ a :=
|
|
begin
|
|
intro Hab,
|
|
have Ha : a, from and.elim_left Hab,
|
|
have Hb : b, from and.elim_right Hab,
|
|
show b ∧ a, from and.intro _ Ha
|
|
end
|