aboutsummaryrefslogtreecommitdiffstats
path: root/examples/switching_input.v
blob: 52261d8f4de453e8ee6c05c06e063ff764979ff7 (plain)
1
2
3
4
5
6
7
8
9
10
Require Import SMTCoq.
Require Import Bool.
Local Open Scope int63_scope.

Parameter m : Z -> Z.
Axiom m_0 : m 0 =? 5.

Lemma cinq_m_0 :
  m 0 =? 5.
Proof. verit_base m_0; vauto. Qed.