Section fsm_experiment.
Inductive state :Type :=
| s1:state
| s2:state.
Inductive input :Type :=
| i1:input
| i2:input.
Definition transitions(s:state)(i:input):state :=
match s, i with
| s1, i1 => s1
| s1, i2 => s2
| s2, i1 => s2
| s2, i2 => s1
end.
Lemma i1_same_state: forall s:state, (transitions s i1) = s.
Proof.
intros.
induction s.
simpl.
reflexivity.
simpl.
reflexivity.
Qed.
Lemma i2_diff_state: forall s:state, (transitions s i2) <> s.
Proof.
intros.
induction s.
simpl.
intuition.
inversion H.
simpl.
intuition.
inversion H.
Qed.
End fsm_experiment.