aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/ideal-features/apply.v
blob: b10d5dbf9c76f0f0737b287e0d2022e16eda28cb (plain)
1
2
3
4
5
6
7
8
9
(* Test propagation of evars from subgoal to brother subgoals *)

(* This does not work (oct 2008) because "match goal" sees "?evar = O" 
   and not "O = O"

Lemma eapply_evar : O=O -> 0=O.
intro H; eapply trans_equal; 
  [apply H | match goal with |- ?x = ?x => reflexivity end].
Qed.