blob: 2d13c0f486fed4099ba0c5bfa0656af95a2d08fd (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
|
(* In order to test the latest thm deps setup, consider this example: *)
theory Depends imports Main begin
lemma I: "A ==> A" and K: "A ==> B ==> A" .
(*
This reports I, K depending on several things; for your internal
dependency graph you may interpret this as each member of {I, K} depending
on all the deps.
*)
end
|