src/HOL/ex/Puzzle.ML
changeset 12486 0ed8bdd883e0
parent 9870 2374ba026fc6
equal deleted inserted replaced
12485:3df60299a6d0 12486:0ed8bdd883e0
    30 Goal "m <= n --> f(m) <= f(n)";
    30 Goal "m <= n --> f(m) <= f(n)";
    31 by (induct_tac "n" 1);
    31 by (induct_tac "n" 1);
    32  by (Simp_tac 1);
    32  by (Simp_tac 1);
    33 by (rtac impI 1);
    33 by (rtac impI 1);
    34 by (etac le_SucE 1);
    34 by (etac le_SucE 1);
    35  by(cut_inst_tac [("n","n")]lemma2 1);
    35  by (cut_inst_tac [("n","n")]lemma2 1);
    36  by(arith_tac 1);
    36  by (arith_tac 1);
    37 by(Asm_simp_tac 1);
    37 by (Asm_simp_tac 1);
    38 qed_spec_mp "f_mono";
    38 qed_spec_mp "f_mono";
    39 
    39 
    40 Goal "f(n) = n";
    40 Goal "f(n) = n";
    41 by (rtac order_antisym 1);
    41 by (rtac order_antisym 1);
    42 by (rtac lemma1 2);
    42 by (rtac lemma1 2);